Issue2756.agda 97 B

1234567891011
  1. module Issue2756 where
  2. module M where
  3. postulate A : Set
  4. module M′ = M
  5. B : Set
  6. B = M′.A