examples.prop_encodableArchive.Examples.PropEncodable

This file has been ported!

Changes since the initial port

The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.

Changes in mathlib3

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(no changes)

(last sync)

Changes in mathlib3port

mathlib3
mathlib3port
Diff
@@ -3,7 +3,7 @@ Copyright (c) 2019 Jeremy Avigad. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Jeremy Avigad
 -/
-import Mathbin.Data.W.Basic
+import Data.W.Basic
 
 #align_import examples.prop_encodable from "leanprover-community/mathlib"@"08b081ea92d80e3a41f899eea36ef6d56e0f1db0"
 
Diff
@@ -2,14 +2,11 @@
 Copyright (c) 2019 Jeremy Avigad. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Jeremy Avigad
-
-! This file was ported from Lean 3 source module examples.prop_encodable
-! leanprover-community/mathlib commit 08b081ea92d80e3a41f899eea36ef6d56e0f1db0
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathbin.Data.W.Basic
 
+#align_import examples.prop_encodable from "leanprover-community/mathlib"@"08b081ea92d80e3a41f899eea36ef6d56e0f1db0"
+
 /-!
 # W types
 
Diff
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Jeremy Avigad
 
 ! This file was ported from Lean 3 source module examples.prop_encodable
-! leanprover-community/mathlib commit 328375597f2c0dd00522d9c2e5a33b6a6128feeb
+! leanprover-community/mathlib commit 08b081ea92d80e3a41f899eea36ef6d56e0f1db0
 ! Please do not edit these lines, except to modify the commit id
 ! if you have ported upstream changes.
 -/
@@ -13,6 +13,9 @@ import Mathbin.Data.W.Basic
 /-!
 # W types
 
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
 The file `data/W.lean` shows that if `α` is an an encodable fintype and for every `a : α`,
 `β a` is encodable, then `W β` is encodable.
 
Diff
@@ -76,16 +76,12 @@ namespace PropForm
 private def constructors (α : Type _) :=
   Sum α (Sum Unit (Sum Unit Unit))
 
--- mathport name: «exprcvar »
 local notation "cvar " a => Sum.inl a
 
--- mathport name: exprcnot
 local notation "cnot" => Sum.inr (Sum.inl Unit.unit)
 
--- mathport name: exprcand
 local notation "cand" => Sum.inr (Sum.inr (Sum.inr Unit.unit))
 
--- mathport name: exprcor
 local notation "cor" => Sum.inr (Sum.inr (Sum.inl Unit.unit))
 
 @[simp]

Changes in mathlib4

mathlib3
mathlib4
style: homogenise porting notes (#11145)

Homogenises porting notes via capitalisation and addition of whitespace.

It makes the following changes:

  • converts "--porting note" into "-- Porting note";
  • converts "porting note" into "Porting note".
Diff
@@ -42,7 +42,7 @@ The next three functions make it easier to construct functions from a small
 `Fin`.
 -/
 
--- porting note: using `![_, _]` notation instead
+-- Porting note: using `![_, _]` notation instead
 #noalign prop_encodable.mk_fn0
 #noalign prop_encodable.mk_fn1
 #noalign prop_encodable.mk_fn2
feat: vertex replacement (#6808)

cliqueFree_of_replaceVertex_cliqueFree is still quite long.

Diff
@@ -30,7 +30,7 @@ show encodability.
 namespace PropEncodable
 
 /-- Propositional formulas with labels from `α`. -/
-inductive PropForm (α : Type _)
+inductive PropForm (α : Type*)
   | var : α → PropForm α
   | not : PropForm α → PropForm α
   | and : PropForm α → PropForm α → PropForm α
@@ -49,7 +49,7 @@ The next three functions make it easier to construct functions from a small
 
 namespace PropForm
 
-private def Constructors (α : Type _) :=
+private def Constructors (α : Type*) :=
   α ⊕ (Unit ⊕ (Unit ⊕ Unit))
 
 local notation "cvar " a => Sum.inl a
@@ -61,13 +61,13 @@ local notation "cand" => Sum.inr (Sum.inr (Sum.inr Unit.unit))
 local notation "cor" => Sum.inr (Sum.inr (Sum.inl Unit.unit))
 
 @[simp]
-private def arity (α : Type _) : Constructors α → Nat
+private def arity (α : Type*) : Constructors α → Nat
   | cvar _ => 0
   | cnot => 1
   | cand => 2
   | cor => 2
 
-variable {α : Type _}
+variable {α : Type*}
 
 instance : ∀ c : Unit ⊕ (Unit ⊕ Unit), NeZero (arity α (.inr c))
   | .inl () => ⟨one_ne_zero⟩
chore: fix grammar mistakes (#6121)
Diff
@@ -11,7 +11,7 @@ import Mathlib.Data.Fin.VecNotation
 /-!
 # W types
 
-The file `Mathlib/Data/W/Basic.lean` shows that if `α` is an an encodable fintype and for every
+The file `Mathlib/Data/W/Basic.lean` shows that if `α` is an encodable fintype and for every
 `a : α`, `β a` is encodable, then `W β` is encodable.
 
 As an example of how this can be used, we show that the type of propositional formulas with
chore: script to replace headers with #align_import statements (#5979)

Open in Gitpod

Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com>

Diff
@@ -2,15 +2,12 @@
 Copyright (c) 2019 Jeremy Avigad. All rights reserved.
 Released under Apache 2.0 license as described in the file LICENSE.
 Authors: Jeremy Avigad
-
-! This file was ported from Lean 3 source module examples.prop_encodable
-! leanprover-community/mathlib commit 328375597f2c0dd00522d9c2e5a33b6a6128feeb
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
 -/
 import Mathlib.Data.W.Basic
 import Mathlib.Data.Fin.VecNotation
 
+#align_import examples.prop_encodable from "leanprover-community/mathlib"@"328375597f2c0dd00522d9c2e5a33b6a6128feeb"
+
 /-!
 # W types
 
chore: tidy various files (#5458)
Diff
@@ -14,8 +14,8 @@ import Mathlib.Data.Fin.VecNotation
 /-!
 # W types
 
-The file `data/W.lean` shows that if `α` is an an encodable fintype and for every `a : α`,
-`β a` is encodable, then `W β` is encodable.
+The file `Mathlib/Data/W/Basic.lean` shows that if `α` is an an encodable fintype and for every
+`a : α`, `β a` is encodable, then `W β` is encodable.
 
 As an example of how this can be used, we show that the type of propositional formulas with
 variables labeled from an encodable type is encodable.
@@ -42,7 +42,7 @@ inductive PropForm (α : Type _)
 
 /-!
 The next three functions make it easier to construct functions from a small
-`fin`.
+`Fin`.
 -/
 
 -- porting note: using `![_, _]` notation instead
chore(Topology/{Paracompact + PartitionOfUnity + Algebra/Order/Compact}): restore a more faithful mathported proof, using the "newer" push_neg (#5132)

These are just three cases where a mathported proof had to be changed, due to unwanted behaviour with push_neg/contradiction. Since #5082 is supposed to fix some issues with these tactics, some of these workarounds can be removed.

Note: this was not in any way systematic, I simply grepped the line after a contra, then grepped for a not and then selected 3 likely candidates. There are potentially more situations like these.

Dependencies 6 + 211

212 files ported (97.2%)
93558 lines ported (97.7%)
Show graph

The unported dependencies are