This repository was archived by the owner on Jul 24, 2024. It is now read-only.
-
Notifications
You must be signed in to change notification settings - Fork 292
[Merged by Bors] - feat(field_theory): finite fields exist #8692
Closed
Closed
Changes from all commits
Commits
Show all changes
40 commits
Select commit
Hold shift + click to select a range
4ee62b2
A first stup
jcommelin c00ee61
char_p
jcommelin b2a56f9
WIP
jcommelin ec29583
adjoin_univ
jcommelin 9b7a8dd
some polynomial lemmas
alexjbest ec8b668
Starting to prove that the first Galois field 'is' zmod p
awainverse 2f45c82
Some more instances, fixed some sorries
awainverse b0556a9
Move one_lt_card
jcommelin d5add51
Some useful lemmas
awainverse 0119513
Merge branch 'finite-fields-exist' of https://github.com/leanprover-c…
awainverse c1a0649
WIP
jcommelin 672a9f7
some refactoring
jcommelin 2513e6a
Merge master.
Ruben-VandeVelde 6ff0478
Fixes
Ruben-VandeVelde 689159e
Attempt proof
Ruben-VandeVelde d20f57a
lemma already in mathlib
alexjbest 9e6c6f6
last sorries?
alexjbest e8c1258
typo
alexjbest 53bd0a5
Fixes
Ruben-VandeVelde 581070c
Apply suggestions from code review
Ruben-VandeVelde 117b6fb
adjust to lemma in mathlib
alexjbest e9fde94
shorter proof
alexjbest b1dedc7
Fix card lemma
Ruben-VandeVelde 8493f99
Merge branch 'finite-fields-exist' of github.com:leanprover-community…
alexjbest d0a11a6
copyright
alexjbest 6d81569
fix names
alexjbest 87c6f30
Move
Ruben-VandeVelde c719b5e
Apply suggestions from code review
Ruben-VandeVelde 10bbba0
Doc
Ruben-VandeVelde 137a6ca
Refactor
Ruben-VandeVelde ce76a53
nicer proof?
alexjbest 3acbe21
Update src/data/zmod/algebra.lean
alexjbest 1744e40
Update algebra.lean
Ruben-VandeVelde 6c5be86
Lint fixes
Ruben-VandeVelde 317527d
Remove card_roots_eq_of_separable_of_splits
Ruben-VandeVelde 8f88967
Move exists_finset_of_splits
Ruben-VandeVelde 0795172
Rename card_eq_pow_finrank
Ruben-VandeVelde a6e03c3
move
Ruben-VandeVelde fdc090d
remove dangerous looking instance
alexjbest de3eef9
oops remove lint
alexjbest File filter
Filter by extension
Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
There are no files selected for viewing
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
| Original file line number | Diff line number | Diff line change |
|---|---|---|
| @@ -0,0 +1,43 @@ | ||
| /- | ||
| Copyright (c) 2021 Johan Commelin. All rights reserved. | ||
| Released under Apache 2.0 license as described in the file LICENSE. | ||
| Authors: Johan Commelin | ||
| -/ | ||
|
|
||
| import data.zmod.basic | ||
| import algebra.algebra.basic | ||
|
|
||
| /-! | ||
| # The `zmod n`-algebra structure on rings whose characteristic divides `n` | ||
| -/ | ||
|
|
||
| namespace zmod | ||
|
|
||
| variables (R : Type*) [ring R] | ||
|
|
||
| section | ||
| variables {n : ℕ} (m : ℕ) [char_p R m] | ||
|
|
||
| /-- The `zmod n`-algebra structure on rings whose characteristic `m` divides `n` -/ | ||
| def algebra' (h : m ∣ n) : algebra (zmod n) R := | ||
| { smul := λ a r, a * r, | ||
| commutes' := λ a r, show (a * r : R) = r * a, | ||
| begin | ||
| rcases zmod.int_cast_surjective a with ⟨k, rfl⟩, | ||
| show zmod.cast_hom h R k * r = r * zmod.cast_hom h R k, | ||
| rw ring_hom.map_int_cast, | ||
| exact commute.cast_int_left r k, | ||
| end, | ||
| smul_def' := λ a r, rfl, | ||
| .. zmod.cast_hom h R } | ||
|
|
||
| end | ||
|
|
||
| section | ||
| variables (n : ℕ) [char_p R n] | ||
|
|
||
| instance : algebra (zmod n) R := algebra' R n (dvd_refl n) | ||
|
|
||
| end | ||
|
|
||
| end zmod | ||
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Oops, something went wrong.
Add this suggestion to a batch that can be applied as a single commit.
This suggestion is invalid because no changes were made to the code.
Suggestions cannot be applied while the pull request is closed.
Suggestions cannot be applied while viewing a subset of changes.
Only one suggestion per line can be applied in a batch.
Add this suggestion to a batch that can be applied as a single commit.
Applying suggestions on deleted lines is not supported.
You must change the existing code in this line in order to create a valid suggestion.
Outdated suggestions cannot be applied.
This suggestion has been applied or marked resolved.
Suggestions cannot be applied from pending reviews.
Suggestions cannot be applied on multi-line comments.
Suggestions cannot be applied while the pull request is queued to merge.
Suggestion cannot be applied right now. Please check back later.
Uh oh!
There was an error while loading. Please reload this page.