Zulip Chat Archive

Stream: general

Topic: recreational group theory


Johan Commelin (May 26 2020 at 06:43):

Exercise A.1.22. The fundamental group of English is generated by the 26 letters a, . . . ,z, subject to all relations w=u where w and u are letter sequences that are pronounced identically in at least some contexts. E.g., gh is trivial since it is silent in some words, and ir = er because of the words “bird” and “her”.

Prove that this group is trivial.

[https://www.math.uni-bielefeld.de/~bux/texts/ggt_notes.pdf]

Mario Carneiro (May 26 2020 at 06:47):

I suppose the goal is to prove that the group is trivial?

Mario Carneiro (May 26 2020 at 06:48):

I wouldn't want to formalize the question though

Johan Commelin (May 26 2020 at 06:50):

No, but you could still prove formally that the group is trivial

Johan Commelin (May 26 2020 at 06:50):

I imagine it would push us towards creating some tools

Mario Carneiro (May 26 2020 at 06:50):

you could prove formally that any group with at least some chosen key subset of relations is trivial

Mario Carneiro (May 26 2020 at 06:50):

but the entire description of the group is quite large

Johan Commelin (May 26 2020 at 06:51):

Well, if we prove that:

G/H is trivial, and H < H', then G/H' is trivial
then I consider that part settled.

Mario Carneiro (May 26 2020 at 06:52):

That still doesn't constitute a formal proof. At the very least you have to write down all the relations and note that the ones you care about are in the list

Mario Carneiro (May 26 2020 at 06:54):

I believe that it is possible to make a convincing argument that there exists in theory a description of a fundamental group of English, and any such description must necessarily contain such and such relations therefore QED, but that's more like a proof of provable statement existence than a proof

Johan Commelin (May 26 2020 at 06:55):

I agree.

Johan Commelin (May 26 2020 at 06:57):

So... the challenge would be: write down an explicit list of relations (like "er" = "ir", with witnesses in the comments), and prove that the free group on 26 letters of the alphabet modulo these relations is trivial.
That is something we can do in principal, but is still nontrivial.

Mario Carneiro (May 26 2020 at 06:57):

that's true

Mario Carneiro (May 26 2020 at 06:58):

I guess I would try to set up the problem such that I need to prove that a = 1, b = 1, ...., z = 1 and conclude

Mario Carneiro (May 26 2020 at 06:58):

with the equalities being regular equalities of elements in a group, so that I can apply cancellation rules as normal

Kevin Buzzard (May 26 2020 at 07:06):

One could also prove the arguably more famous theorem of Zagier at al, where two words are the same if they're pronounced the same way. They proved that the homophonic group was trivial for English and French IIRC

Kevin Buzzard (May 26 2020 at 07:07):

https://projecteuclid.org/euclid.em/1062620828

Kevin Buzzard (May 26 2020 at 07:08):

This is the same journal that will have a maths formalisation issue next year

Scott Morrison (May 26 2020 at 07:15):

"One could give a proof with a more topological flavor of the triviality of f using cerf = serre."

Kevin Buzzard (May 26 2020 at 07:17):

I remember this caused quite a stir when it came out

Mario Carneiro (May 26 2020 at 07:35):

huh, there seem to be a lot of missing theorems here around free_group and presented_group

Mario Carneiro (May 26 2020 at 07:36):

it isn't even proven that the relations in a presented group are trivialized in the group

Mario Carneiro (May 26 2020 at 07:36):

also universal properties in terms of membership in a subgroup

Kevin Buzzard (May 26 2020 at 07:53):

I think formalising this theorem would (a) be easy (b) be interesting and (c) teach us about holes in mathlib

Kevin Buzzard (May 26 2020 at 07:54):

It would probably also be something which undergraduates could do and send to Exp Math :-)

Mario Carneiro (May 26 2020 at 07:59):

import group_theory.presented_group

namespace free_group

theorem subgroup_induction {α} {p : set (free_group α)} [is_subgroup p]
  (h :  a, of a  p) (x : free_group α) : x  p :=
free_group.induction_on x is_submonoid.one_mem h
  (λ _, is_subgroup.inv_mem) (λ _ _, is_submonoid.mul_mem)

end free_group

namespace english

inductive alphabet
| a | b | c | d | e | f | g | h | i | j | k | l | m
| n | o | p | q | r | s | t | u | v | w | x | y | z

section
open alphabet
open free_group (of)

inductive rel : free_group alphabet  free_group alphabet  Prop
| er_ir : rel (of e * of r) (of i * of r)
| gh_ : rel (of g * of h) 1
-- add relations here
end

@[derive group]
def G := presented_group {z |  x y, rel x y  z = x⁻¹ * y}
instance : has_coe alphabet G := presented_group.of

theorem to_G {a b : free_group alphabet} (h : rel a b) :
  (quotient_group.mk a : G) = quotient_group.mk b :=
quotient_group.eq.2 (group.subset_normal_closure a, b, h, rfl)

open alphabet
theorem foo (γ : G) : γ = 1 :=
begin
  suffices :  α : alphabet, (α : G) = 1,
  { refine quotient_group.induction_on' γ (λ z, _),
    refine (@is_group_hom.mem_ker _ _ _ quotient_group.mk z).1 _,
    refine free_group.subgroup_induction _ z,
    intro, rw is_group_hom.mem_ker, exact this _ },
  clear γ, intro α,
  have : (e * r : G) = i * r := to_G rel.er_ir,
  have : (g * h : G) = 1 := to_G rel.gh_,
  cases α,
  -- have fun
end

end english

Kenny Lau (May 26 2020 at 09:44):

Kenny Lau (May 26 2020 at 09:45):

til "halfpenny" is pronounced /ˈheɪp(ə)ni/ ???

Mario Carneiro (May 26 2020 at 09:45):

ha-penny

Sebastien Gouezel (May 26 2020 at 09:46):

What is fivepence, and how is it pronounced?

Mario Carneiro (May 26 2020 at 09:46):

fi-pence I think

Kenny Lau (May 26 2020 at 09:46):

@Kevin Buzzard please fix your language

Sebastien Gouezel (May 26 2020 at 09:46):

Come on, they are even more crazy than I thought.

Mario Carneiro (May 26 2020 at 09:46):

I question the monsieur example though

Mario Carneiro (May 26 2020 at 09:47):

I get something like n = õ - o

Kenny Lau (May 26 2020 at 09:47):

how about "hymn"

Kenny Lau (May 26 2020 at 09:47):

there's no nasalization in "monsieur" though

Kenny Lau (May 26 2020 at 09:48):

not even in French

Chris Hughes (May 26 2020 at 09:48):

aar=araar = ar because of aardvark and car, so a=1a = 1
mb=mmb = m because of plumb and plum so b=1b = 1
ck=kck = k because of back and book so c=1c = 1
d=1d = 1
ea=aea = a because of bread and bed so e=1e = 1
f=1f = 1 because of Ffion and Fiona
g=1g = 1 because it is silent in Gnasher
h=1h = 1 because it is silent in hour
i=eei = ee because of ski and bee, so i=1i=1
j=1j=1 because g=1g=1 and page and Japan
$$k = 1$ since it is silent in knife
l=1l=1 because of nil and
m=1m=1 because it is silent in mnemonic
n=1n=1 because it is silent in autumn
oo=ooo = o because of tomb and boom
p=1p=1 because it is silent in pneumatic
q=cq = c because of quarter and cat, so q=1q=1
ar=aar = a because of grass and car so r=1r = 1 (South East England specific)
s=cs=c because of ceiling, so s=1s=1
t=1t=1 because it is silent in castle
u=oou=oo because of flu and boo sso u=1u=1
v=1v=1
ow=oeow=oe because of tow and toe, so w=1w=1
x=cksx = cks because of fox and kicks, so x=1x = 1
y=eey=ee because of quickly and bee, so y=1y=1
z=xz = x because of xylophone so z=1z=1

Kenny Lau (May 26 2020 at 09:48):

@Sebastien Gouezel can confirm

Chris Hughes (May 26 2020 at 09:48):

I was stuck on dd and vv

Patrick Massot (May 26 2020 at 09:48):

The French pronunciation of monsieur is completely random, as often happen with very common words (they are used a lot, hence in bad shape)

Johan Commelin (May 26 2020 at 09:49):

Is rijsttafel an English word?

Patrick Massot (May 26 2020 at 09:49):

sounds like Dutch to me

Mario Carneiro (May 26 2020 at 09:49):

aha, as in it sounds like "misier"

Mario Carneiro (May 26 2020 at 09:49):

it is definitely dutch

Mario Carneiro (May 26 2020 at 09:50):

well, it's a dutch word for an indonesian meal

Chris Hughes (May 26 2020 at 09:50):

fivepence is cheating. There must be a better one for vv

Kenny Lau (May 26 2020 at 09:50):

revving?

Kenny Lau (May 26 2020 at 09:50):

for d how about add

Chris Hughes (May 26 2020 at 09:51):

I feel like double letters in the middle of words makes it too easy.

Kenny Lau (May 26 2020 at 09:52):

all vowels are equivalent because they all get reduced

Sebastien Gouezel (May 26 2020 at 09:52):

Chris Hughes said:

p=1p=1 because it is silent in pneumatic

What?

Kenny Lau (May 26 2020 at 09:53):

yeah it's also silent in pterodactyl

Kenny Lau (May 26 2020 at 09:53):

and psychology

Kevin Buzzard (May 26 2020 at 09:53):

I have never heard of the word fivepence and have no idea about this missing v

Sebastien Gouezel (May 26 2020 at 09:54):

I knew about psychology, I guess the other ones are less common.

Kenny Lau (May 26 2020 at 09:54):

how are you supposed to pronounce "pn" in french

Kevin Buzzard (May 26 2020 at 09:54):

But "hay-p'ny" for halfpenny was common when that coin existed (it disappeared in the mid 80s)

Kenny Lau (May 26 2020 at 09:55):

D is shirking its auditory duties in handkerchief and mostly doing the same in handsome. Its appearance in Wednesday can only be seen as some kind of cruel joke.

Patrick Massot (May 26 2020 at 09:55):

In French pneumatique uses both the p and n

Kenny Lau (May 26 2020 at 09:55):

is "Wednesday" cheating?

Kenny Lau (May 26 2020 at 09:55):

how about "Godmanchester" (pronounced "Gumster")

Patrick Massot (May 26 2020 at 09:56):

Wednesday seems totally fair

Kenny Lau (May 26 2020 at 09:56):

there's a silent d, silent n, silent ch

Chris Hughes (May 26 2020 at 09:56):

I knew someone who lived in Godmanchester and he didn't say Gumster

Patrick Massot (May 26 2020 at 09:56):

City names are cheating

Kenny Lau (May 26 2020 at 09:57):

V is at this point the only letter that refuses to be unheard in any established word of the language. And yet a dark cloud gathers on the horizon: in late May 2017 a much-followed and likely sleep-addled Twitter user tweeted out what was clearly a partially developed composition. The Internet seized on the enigmatic final word and discussed it ad nauseam. Of the myriad pronunciations suggested for this non-word, several of the strongest contenders had a silent v.

Kenny Lau (May 26 2020 at 09:57):

so Merriam Webster doesn't have any better for v

Kenny Lau (May 26 2020 at 09:57):

that just means it can't be silent

Kenny Lau (May 26 2020 at 09:57):

it can still be related via non-trivial means

Chris Hughes (May 26 2020 at 09:58):

But I can't think of words where any other letter is pronounced vv either.

Kenny Lau (May 26 2020 at 09:58):

I feel like the closest would be some German borrowings where the "v" is pronounced "f"

Amelia Livingston (May 26 2020 at 10:00):

of?

Kenny Lau (May 26 2020 at 10:00):

Some of you may be happy to know that we have at this point only one English word in which the j is silent: marijuana.

Kenny Lau (May 26 2020 at 10:04):

@Chris Hughes your example for e is invalid: it only shows ea=e, i.e. a=1

Chris Hughes (May 26 2020 at 10:05):

Oops.

Kenny Lau (May 26 2020 at 10:05):

how about meat = meet

Chris Hughes (May 26 2020 at 10:05):

That works.

Chris Hughes (May 26 2020 at 10:05):

Maybe a better example for F would be good as well.

Kenny Lau (May 26 2020 at 10:06):

and for f how about cough

Rob Lewis (May 26 2020 at 10:07):

Mario Carneiro said:

well, it's a dutch word for an indonesian meal

It's a Dutch word for Indonesian food served in a style unique to the Netherlands, or at least I've been told. You all ate this at Lean Together 2019 ;)

Kenny Lau (May 26 2020 at 10:20):

(largely based on Chris' answer)
a: bread / bred
b: plumb
c: scene / seen
d: Wednesday
e: meat / meet
f: cough
g: gnash
h: hour
i: business
j: Japan / page
k: knife
l: salmon
m: mnemonic
n: autumn
o: people
p: psychology
q: pique / peek
r: forecastle (pronounced "foe-ksel"???)
s: seed / cede
t: listen
u: guard
v: of
w: write / rite
x: xylophone (z)
y: sky / tie
z: disaster (s)

Chris Hughes (May 26 2020 at 10:25):

Never heard of forecastle

Kenny Lau (May 26 2020 at 10:27):

The forecastle (/ˈfoʊksəl/ FOHK-səl; abbreviated fo'c'sle or fo'c's'le) is the upper deck of a sailing ship forward of the foremast, or the forward part of a ship with the sailors' living quarters.

Chris Hughes (May 26 2020 at 10:28):

That'll be why I haven't heard of it. I'm not an 18th century sailor.

Patrick Stevens (May 26 2020 at 12:17):

In a similar vein you can get "rollock" and "rowlock" which are pronounced the same way

Patrick Stevens (May 26 2020 at 12:17):

Lots of good nautical words


Last updated: Dec 20 2023 at 11:08 UTC