@@ -192,11 +192,11 @@ private
192192 ⊤ ∧ y ≈⟨ ∧-identityˡ _ ⟩
193193 y ∎
194194
195- ⊥≉ ⊤ : ¬ ⊥ ≈ ⊤
196- ⊥≉ ⊤ = lemma ⊥ ⊤ (∧-identityʳ _) (∨-zeroʳ _)
195+ ¬⊥≈ ⊤ : ¬ ⊥ ≈ ⊤
196+ ¬⊥≈ ⊤ = lemma ⊥ ⊤ (∧-identityʳ _) (∨-zeroʳ _)
197197
198- ⊤≉ ⊥ : ¬ ⊤ ≈ ⊥
199- ⊤≉ ⊥ = lemma ⊤ ⊥ (∧-zeroʳ _) (∨-identityʳ _)
198+ ¬⊤≈ ⊥ : ¬ ⊤ ≈ ⊥
199+ ¬⊤≈ ⊥ = lemma ⊤ ⊥ (∧-zeroʳ _) (∨-identityʳ _)
200200
201201¬-involutive : Involutive ¬_
202202¬-involutive x = lemma (¬ x) x (∧-complementˡ _) (∨-complementˡ _)
@@ -308,7 +308,7 @@ module XorRing
308308 ⊕-identityˡ x = begin
309309 ⊥ ⊕ x ≈⟨ ⊕-def _ _ ⟩
310310 (⊥ ∨ x) ∧ ¬ (⊥ ∧ x) ≈⟨ helper (∨-identityˡ _) (∧-zeroˡ _) ⟩
311- x ∧ ¬ ⊥ ≈⟨ ∧-congˡ ⊥≉ ⊤ ⟩
311+ x ∧ ¬ ⊥ ≈⟨ ∧-congˡ ¬⊥≈ ⊤ ⟩
312312 x ∧ ⊤ ≈⟨ ∧-identityʳ _ ⟩
313313 x ∎
314314
@@ -536,3 +536,23 @@ _⊕_ : Op₂ Carrier
536536x ⊕ y = (x ∨ y) ∧ ¬ (x ∧ y)
537537
538538module DefaultXorRing = XorRing _⊕_ (λ _ _ → refl)
539+
540+
541+ ------------------------------------------------------------------------
542+ -- DEPRECATED NAMES
543+ ------------------------------------------------------------------------
544+ -- Please use the new names as continuing support for the old names is
545+ -- not guaranteed.
546+
547+ -- Version 2.3
548+
549+ ⊥≉⊤ = ¬⊥≈⊤
550+ {-# WARNING_ON_USAGE ⊥≉⊤
551+ "Warning: ⊥≉⊤ was deprecated in v2.3.
552+ Please use ¬⊥≈⊤ instead."
553+ #-}
554+ ⊤≉⊥ = ¬⊤≈⊥
555+ {-# WARNING_ON_USAGE ⊤≉⊥
556+ "Warning: ⊤≉⊥ was deprecated in v2.3.
557+ Please use ¬⊤≈⊥ instead."
558+ #-}
0 commit comments