File tree Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -297,8 +297,8 @@ record Semigroup : Set (suc (a ⊔ ℓ)) where
297297-- laws. These correspond more or less to what the definitions would
298298-- be in non-dependently typed languages like Haskell.
299299
300- -- Each bundle thereofre has a corresponding raw bundle that only
301- -- include the laws but not the operations .
300+ -- Each bundle therefore has a corresponding raw bundle that only
301+ -- includes the operations, but not the laws .
302302
303303record RawMagma c ℓ : Set (suc (c ⊔ ℓ)) where
304304 infixl 7 _∙_
@@ -328,9 +328,9 @@ record RawMonoid c ℓ : Set (suc (c ⊔ ℓ)) where
328328total⇒refl : ∀ {_∼_ : Rel A ℓ} → Total _∼_ → Reflexive _∼_
329329total⇒refl = {!!}
330330
331- idˡ+ comm⇒idʳ : ∀ {_≈_ : Rel A ℓ} {e _∙_} → Commutative _≈_ _∙_ →
331+ idˡ∧ comm⇒idʳ : ∀ {_≈_ : Rel A ℓ} {e _∙_} → Commutative _≈_ _∙_ →
332332 LeftIdentity _≈_ e _∙_ → RightIdentity _≈_ e _∙_
333- idˡ+ comm⇒idʳ = {!!}
333+ idˡ∧ comm⇒idʳ = {!!}
334334
335335------------------------------------------------------------------------
336336-- X.Construct
You can’t perform that action at this time.
0 commit comments